src/HOL/ex/Tree23.thy
changeset 55414 eab03e9cee8a
parent 55413 a8e96847523c
child 55417 01fbfb60c33e
equal deleted inserted replaced
55413:a8e96847523c 55414:eab03e9cee8a
   330 "dfull n (Some (p, (False, t'))) \<longleftrightarrow> full (Suc n) t'"
   330 "dfull n (Some (p, (False, t'))) \<longleftrightarrow> full (Suc n) t'"
   331 
   331 
   332 lemmas dfull_case_intros =
   332 lemmas dfull_case_intros =
   333   ord.exhaust [where y=y and P="dfull a (ord_case b c d y)"]
   333   ord.exhaust [where y=y and P="dfull a (ord_case b c d y)"]
   334   option.exhaust [of y "dfull a (case_option b c y)"]
   334   option.exhaust [of y "dfull a (case_option b c y)"]
   335   prod.exhaust [where y=y and P="dfull a (prod_case b y)"]
   335   prod.exhaust [of y "dfull a (case_prod b y)"]
   336   bool.exhaust [where y=y and P="dfull a (bool_case b c y)"]
   336   bool.exhaust [of y "dfull a (case_bool b c y)"]
   337   tree23.exhaust [where y=y and P="dfull a (Some (b, tree23_case c d e y))"]
   337   tree23.exhaust [where y=y and P="dfull a (Some (b, tree23_case c d e y))"]
   338   tree23.exhaust [where y=y and P="full a (tree23_case b c d y)"]
   338   tree23.exhaust [where y=y and P="full a (tree23_case b c d y)"]
   339   for a b c d e y
   339   for a b c d e y
   340 
   340 
   341 lemma dfull_del: "full (Suc n) t \<Longrightarrow> dfull n (del k t)"
   341 lemma dfull_del: "full (Suc n) t \<Longrightarrow> dfull n (del k t)"