src/HOL/ex/Multiquote.thy
changeset 8627 44ec33bb5c5b
parent 8578 3b9e3c782eb2
child 9297 bafe45732b10
equal deleted inserted replaced
8626:76e3913ff421 8627:44ec33bb5c5b
    38 
    38 
    39 text {* advanced examples *};
    39 text {* advanced examples *};
    40 term ".(.(` `x + `y).).";
    40 term ".(.(` `x + `y).).";
    41 term ".(.(` `x + `y). o `f).";
    41 term ".(.(` `x + `y). o `f).";
    42 term ".(`(f o `g)).";
    42 term ".(`(f o `g)).";
    43 term ".(.(`(`(f o `g))).).";
    43 term ".(.( ` `(f o `g) ).).";
    44 
    44 
    45 end;
    45 end;