Quot/Examples/AbsRepTest.thy
changeset 922 a2589b4bc442
parent 918 7be9b054f672
child 1097 551eacf071d7
equal deleted inserted replaced
921:dae038c8cd69 922:a2589b4bc442
     1 theory AbsRepTest
     1 theory AbsRepTest
     2 imports "../QuotMain" "../QuotList" "../QuotOption" "../QuotSum" "../QuotProd" List
     2 imports "../QuotMain" "../QuotList" "../QuotOption" "../QuotSum" "../QuotProd" List
     3 begin
     3 begin
     4 
     4 
       
     5 
       
     6 (*
     5 ML_command "ProofContext.debug := false"
     7 ML_command "ProofContext.debug := false"
     6 ML_command "ProofContext.verbose := false"
     8 ML_command "ProofContext.verbose := false"
       
     9 *)
     7 
    10 
     8 ML {*
    11 ML {*
     9 val ctxt0 = @{context}
    12 val ctxt0 = @{context}
    10 val ty = Syntax.read_typ ctxt0 "bool"  
    13 val ty = Syntax.read_typ ctxt0 "bool"  
    11 val ctxt1 = Variable.declare_typ ty ctxt0 
    14 val ctxt1 = Variable.declare_typ ty ctxt0