src/HOL/BNF/Ctr_Sugar.thy
changeset 56013 d64a4ef26edb
parent 56012 cfb21e03fe2a
parent 56008 30666a281ae3
child 56014 748778ac0ab8
     1.1 --- a/src/HOL/BNF/Ctr_Sugar.thy	Thu Dec 05 17:52:12 2013 +0100
     1.2 +++ /dev/null	Thu Jan 01 00:00:00 1970 +0000
     1.3 @@ -1,30 +0,0 @@
     1.4 -(*  Title:      HOL/BNF/Ctr_Sugar.thy
     1.5 -    Author:     Jasmin Blanchette, TU Muenchen
     1.6 -    Copyright   2012
     1.7 -
     1.8 -Wrapping existing freely generated type's constructors.
     1.9 -*)
    1.10 -
    1.11 -header {* Wrapping Existing Freely Generated Type's Constructors *}
    1.12 -
    1.13 -theory Ctr_Sugar
    1.14 -imports Main
    1.15 -keywords
    1.16 -  "wrap_free_constructors" :: thy_goal and
    1.17 -  "no_discs_sels" and
    1.18 -  "rep_compat"
    1.19 -begin
    1.20 -
    1.21 -lemma iffI_np: "\<lbrakk>x \<Longrightarrow> \<not> y; \<not> x \<Longrightarrow> y\<rbrakk> \<Longrightarrow> \<not> x \<longleftrightarrow> y"
    1.22 -by (erule iffI) (erule contrapos_pn)
    1.23 -
    1.24 -lemma iff_contradict:
    1.25 -"\<not> P \<Longrightarrow> P \<longleftrightarrow> Q \<Longrightarrow> Q \<Longrightarrow> R"
    1.26 -"\<not> Q \<Longrightarrow> P \<longleftrightarrow> Q \<Longrightarrow> P \<Longrightarrow> R"
    1.27 -by blast+
    1.28 -
    1.29 -ML_file "Tools/ctr_sugar_util.ML"
    1.30 -ML_file "Tools/ctr_sugar_tactics.ML"
    1.31 -ML_file "Tools/ctr_sugar.ML"
    1.32 -
    1.33 -end