Theory Pairing_Heap_Tree_Analysis2

(* Author: Hauke Brinkop and Tobias Nipkow *)

section ‹Pairing Heaps›

subsection ‹Binary Tree Representation›

theory Pairing_Heap_Tree_Analysis2
imports  
  Pairing_Heap.Pairing_Heap_Tree
  Amortized_Framework
  Priority_Queue_ops_merge
  Lemmas_log
begin

text
‹Verification of logarithmic bounds on the amortized complexity of pairing heaps.
As in cite"FredmanSST86" and "Brinkop", except that the treatment of @{const pass1} is simplified.
TODO: convert the other Pairing Heap analyses to this one.›

fun len :: "'a tree  nat" where 
  "len Leaf = 0"
| "len (Node _ _ r) = 1 + len r"

fun Φ :: "'a tree  real" where
  "Φ Leaf = 0"
| "Φ (Node l x r) = log 2 (size (Node l x r)) + Φ l + Φ r"

lemma link_size[simp]: "size (link hp) = size hp" 
  by (cases hp rule: link.cases) simp_all

lemma size_pass1: "size (pass1 hp) = size hp" 
  by (induct hp rule: pass1.induct) simp_all

lemma size_pass2: "size (pass2 hp) = size hp" 
  by (induct hp rule: pass2.induct) simp_all

lemma size_merge: 
  "is_root h1  is_root h2  size (merge h1 h2) = size h1 + size h2"
  by (simp split: tree.splits)

lemma ΔΦ_insert: "is_root hp  Φ (insert x hp) - Φ hp  log 2  (size hp + 1)"
  by (simp split: tree.splits)

lemma ΔΦ_merge:
  assumes "h1 = Node hs1 x1 Leaf" "h2 = Node hs2 x2 Leaf" 
  shows "Φ (merge h1 h2) - Φ h1 - Φ h2  log 2 (size h1 + size h2) + 1" 
proof -
  let ?hs = "Node hs1 x1 (Node hs2 x2 Leaf)"
  have "Φ (merge h1 h2) = Φ (link ?hs)" using assms by simp
  also have " = Φ hs1 + Φ hs2 + log 2 (size hs1 + size hs2 + 1) + log 2 (size hs1 + size hs2 + 2)"
    by (simp add: algebra_simps)
  also have " = Φ hs1 + Φ hs2 + log 2 (size hs1 + size hs2 + 1) + log 2 (size h1 + size h2)"
     using assms by simp
  finally have "Φ (merge h1 h2) = " .
  have "Φ (merge h1 h2) - Φ h1 - Φ h2 =
   log 2 (size hs1 + size hs2 + 1) + log 2 (size h1 + size h2)
   - log 2 (size hs1 + 1) - log 2 (size hs2 + 1)"
     using assms by (simp add: algebra_simps)
  also have "  log 2 (size h1 + size h2) + 1"
    using ld_le_2ld[of "size hs1" "size hs2"] assms by (simp add: algebra_simps)
  finally show ?thesis .
qed

lemma ΔΦ_pass1: "Φ (pass1 hs) - Φ hs   2 * log 2 (size hs + 1) - len hs + 2"
proof (induction hs rule: pass1.induct)
  case (1 hs1 x hs2 y hs)
  let ?h = "Node hs1 x (Node hs2 y hs)"
  let ?n1 = "size hs1"
  let ?n2 = "size hs2" let ?m = "size hs"
  have "Φ (pass1 ?h) - Φ ?h = Φ (pass1 hs) + log 2 (?n1+?n2+1) - Φ hs - log 2 (?n2+?m+1)" 
    by (simp add: size_pass1 algebra_simps)
  also have "  log 2 (?n1+?n2+1) - log 2 (?n2+?m+1) + 2 * log 2 (?m + 1) - len hs + 2" 
    using "1.IH" by (simp)
  also have "  2 * log 2 (?n1+?n2+?m+2) - log 2 (?n2+?m+1) + log 2 (?m + 1) - len hs" 
        using ld_sum_inequality [of "?n1+?n2+1" "?m + 1"] by(simp)
  also have "  2 * log 2 (?n1+?n2+?m+2) - len hs" by simp
  also have " = 2 * log 2 (size ?h) - len ?h + 2" by simp
  also have "  2 * log 2 (size ?h + 1) - len ?h + 2" by simp
  finally show ?case .
qed simp_all

lemma ΔΦ_pass2: "hs  Leaf  Φ (pass2 hs) - Φ hs  log 2 (size hs)"
proof (induction hs)
  case (Node hs1 x hs)
  thus ?case 
  proof (cases hs)
    case 1: (Node hs2 y r)
    let ?h = "Node hs1 x hs"
    obtain hs3 a where 2: "pass2 hs = Node hs3 a Leaf" 
      using pass2_struct 1 by force
    hence 3: "size hs = size " using size_pass2 by metis
    have link: "Φ(link(Node hs1 x (pass2 hs))) - Φ hs1 - Φ (pass2 hs) =
          log 2 (size hs1 + size hs + 1) + log 2 (size hs1 + size hs) - log 2 (size hs)"
      using 2 3 by (simp add: algebra_simps)
    have "Φ (pass2 ?h) - Φ ?h =
        Φ (link (Node hs1 x (pass2 hs))) - Φ hs1 - Φ hs - log 2 (size hs1 + size hs + 1)"
      by (simp)
    also have " = Φ (pass2 hs) - Φ hs + log 2 (size hs1 + size hs) - log 2 (size hs)"
      using link by linarith
    also have "  log 2 (size hs1 + size hs)"
      using Node.IH(2) 1 by simp
    also have "  log 2 (size ?h)" using 1 by simp
    finally show ?thesis .
  qed simp
qed simp

corollary ΔΦ_pass2': "Φ (pass2 hs) - Φ hs  log 2 (size hs + 1)"
proof cases
  assume "hs = Leaf" thus ?thesis by simp
next
  assume "hs  Leaf"
  hence "log 2 (size hs)  log 2 (size hs + 1)" using eq_size_0 by fastforce
  then show ?thesis using ΔΦ_pass2[OF hs  Leaf] by linarith
qed

lemma ΔΦ_del_min:
  "Φ (del_min (Node hs x Leaf)) - Φ (Node hs x Leaf) 
   2 * log 2 (size hs + 1) - len hs + 2"
proof -
  have "Φ (del_min (Node hs x Leaf)) - Φ (Node hs x Leaf) =
        Φ (pass2 (pass1 hs)) - (log 2 (1 + real (size hs)) + Φ hs)" by simp
  also have "  Φ (pass1 hs) - Φ hs"
    using ΔΦ_pass2' [of "pass1 hs"] by(simp add: size_pass1)
  also have "  2 * log 2 (size hs + 1) - len hs + 2" by(rule ΔΦ_pass1)
  finally show ?thesis .
qed

lemma is_root_merge:
  "is_root h1  is_root h2  is_root (merge h1 h2)"
by (simp split: tree.splits)

lemma is_root_insert: "is_root h  is_root (insert x h)"
by (simp split: tree.splits)

lemma is_root_del_min:
  assumes "is_root h" shows "is_root (del_min h)"
proof (cases h)
  case [simp]: (Node hs1 x hs)
  have "hs = Leaf" using assms by simp
  thus ?thesis 
  proof (cases hs1)
    case (Node hs2 y hs')
    then obtain la a ra where "pass1 hs1 = Node a la ra" 
      using pass1_struct by blast
    moreover obtain lb b where "pass2  = Node b lb Leaf"
      using pass2_struct by blast
    ultimately show ?thesis using assms by simp
  qed simp
qed simp

lemma pass1_len: "len (pass1 h)  len h"
by (induct h rule: pass1.induct) simp_all

fun exec :: "'a :: linorder op  'a tree list  'a tree" where
"exec Empty [] = Leaf" | 
"exec Del_min [h] = del_min h" |
"exec (Insert x) [h] = insert x h" |
"exec Merge [h1,h2] = merge h1 h2"

fun T_pass1 :: "'a tree  nat" where
"T_pass1 (Node _ _ (Node _ _ hs')) = T_pass1 hs' + 1" |
"T_pass1 h = 1"

fun T_pass2 :: "'a tree  nat" where
  "T_pass2 Leaf = 1"
| "T_pass2 (Node _ _ hs) = T_pass2 hs + 1"

fun T_del_min :: "('a::linorder) tree  nat" where
"T_del_min Leaf = 1" |
"T_del_min (Node hs _ _) = T_pass2 (pass1 hs) + T_pass1 hs + 1"

fun T_insert :: "'a  'a tree  nat" where
"T_insert a h = 1"

fun T_merge :: "'a tree  'a tree  nat" where
"T_merge h1 h2 = 1"

lemma A_del_min: assumes "is_root h"
shows "T_del_min h + Φ(del_min h) - Φ h  2 * log 2 (size h + 1) + 5"
proof (cases h)
  case [simp]: (Node hs1 x hs)
  have "T_pass2 (pass1 hs1) + real(T_pass1 hs1)  real(len hs1) + 2"
    by (induct hs1 rule: pass1.induct) simp_all
  moreover have "Φ (del_min h) - Φ h  2 * log 2 (size h + 1) - len hs1 + 2"
  proof -
    have "Φ (del_min h) - Φ h  2 * log 2 (size hs1 + 1) - len hs1 + 2"
      using  ΔΦ_del_min[of "hs1" "x"] assms by simp
    also have "  2 * log 2 (size h + 1) - len hs1 + 2" by fastforce
    finally show ?thesis .
  qed
  ultimately show ?thesis by(simp)
qed simp

lemma A_insert: "is_root h  T_insert a h + Φ(insert a h) - Φ h  log 2 (size h + 1) + 1"
by(drule ΔΦ_insert) simp

lemma A_merge: assumes "is_root h1" "is_root h2"
shows "T_merge h1 h2 + Φ(merge h1 h2) - Φ h1 - Φ h2  log 2 (size h1 + size h2 + 1) + 2"
proof (cases h1)
  case Leaf thus ?thesis by (cases h2) auto
next
  case h1: Node
  show ?thesis
  proof (cases h2)
    case Leaf thus ?thesis using h1 by simp
  next
    case h2: Node
    have "Φ (merge h1 h2) - Φ h1 - Φ h2  log 2 (real (size h1 + size h2)) + 1"
      apply(rule ΔΦ_merge) using h1 h2 assms by auto
    also have "  log 2 (size h1 + size h2 + 1) + 1" by (simp add: h1)
    finally show ?thesis by(simp add: algebra_simps)
  qed
qed

fun cost :: "'a :: linorder op  'a tree list  nat" where
  "cost Empty [] = 1"
| "cost Del_min [h] = T_del_min h"
| "cost (Insert a) [h] = T_insert a h"
| "cost Merge [h1,h2] = T_merge h1 h2"

fun U :: "'a :: linorder op  'a tree list  real" where
  "U Empty [] = 1"
| "U (Insert a) [h] = log 2 (size h + 1) + 1"
| "U Del_min [h] = 2 * log 2 (size h + 1) + 5"
| "U Merge [h1,h2] = log 2 (size h1 + size h2 + 1) + 2"

interpretation Amortized
where arity = arity and exec = exec and cost = cost and inv = is_root 
and Φ = Φ and U = U
proof (standard, goal_cases)
  case (1 _ f) thus ?case using is_root_insert is_root_del_min is_root_merge
    by (cases f) (auto simp: numeral_eq_Suc)
next
  case (2 s) show ?case by (induct s) simp_all
next
  case (3 ss f) show ?case 
  proof (cases f)
    case Empty with 3 show ?thesis by(auto)
  next
    case Insert
    then obtain h where "ss = [h]" "is_root h" using 3 by auto
    thus ?thesis using Insert ΔΦ_insert 3 by auto
  next
    case Del_min
    then obtain h where [simp]: "ss = [h]" using 3 by auto
    show ?thesis using A_del_min[of h] 3 Del_min by simp
  next
    case Merge
    then obtain h1 h2 where "ss = [h1,h2]" "is_root h1" "is_root h2"
      using 3 by (auto simp: numeral_eq_Suc)
    with A_merge[of h1 h2] Merge show ?thesis by simp
  qed
qed

end