src/Doc/Tutorial/Types/Axioms.thy
changeset 72991 d0a0b74f0ad7
parent 69597 ff784d5a5bfb
child 76987 4c275405faae
equal deleted inserted replaced
72990:db8f94656024 72991:d0a0b74f0ad7
     1 (*<*)theory Axioms imports Overloading Setup begin(*>*)
     1 (*<*)theory Axioms imports Overloading "../Setup" begin(*>*)
     2 
     2 
     3 subsection \<open>Axioms\<close>
     3 subsection \<open>Axioms\<close>
     4 
     4 
     5 text \<open>Attaching axioms to our classes lets us reason on the level of
     5 text \<open>Attaching axioms to our classes lets us reason on the level of
     6 classes.  The results will be applicable to all types in a class, just
     6 classes.  The results will be applicable to all types in a class, just