1.1 --- a/src/HOL/Extraction.thy Mon Apr 06 22:11:01 2015 +0200
1.2 +++ b/src/HOL/Extraction.thy Mon Apr 06 23:14:05 2015 +0200
1.3 @@ -34,8 +34,8 @@
1.4 True_implies_equals TrueE
1.5
1.6 lemmas [extraction_expand_def] =
1.7 - induct_forall_def induct_implies_def induct_equal_def induct_conj_def
1.8 - induct_true_def induct_false_def
1.9 + HOL.induct_forall_def HOL.induct_implies_def HOL.induct_equal_def HOL.induct_conj_def
1.10 + HOL.induct_true_def HOL.induct_false_def
1.11
1.12 datatype (plugins only: code extraction) sumbool = Left | Right
1.13